c50227ea6e
This commit also adds the tactic rapply that corresponds to the previous semantics we have been using.
14 lines
376 B
Text
14 lines
376 B
Text
import logic
|
|
open bool eq.ops tactic
|
|
|
|
constants a b c : bool
|
|
axiom H1 : a = b
|
|
axiom H2 : b = c
|
|
|
|
check show a = c, from H1 ⬝ H2
|
|
print "------------"
|
|
check have e1 [visible] : a = b, from H1,
|
|
have e2 : a = c, by apply eq.trans; apply e1; apply H2,
|
|
have e3 : c = a, from e2⁻¹,
|
|
have e4 [visible] : b = a, from e1⁻¹,
|
|
show b = c, from e1⁻¹ ⬝ e2
|