cbc81ea6c5
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
9 lines
249 B
Text
9 lines
249 B
Text
import logic
|
|
using tactic
|
|
|
|
definition my_tac := repeat ([ apply @and_intro
|
|
| apply @refl
|
|
])
|
|
tactic_hint my_tac
|
|
|
|
theorem T1 {A : Type} {B : Type} (a : A) (b c : B) : a = a ∧ b = b ∧ c = c
|