4946f55290
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
21 lines
339 B
Text
21 lines
339 B
Text
import logic
|
|
open eq
|
|
section
|
|
parameter {A : Type}
|
|
theorem T {a b : A} (H : a = b) : b = a
|
|
:= symm H
|
|
parameters x y : A
|
|
hypothesis H : x = y
|
|
check T H
|
|
check T
|
|
end
|
|
|
|
section
|
|
parameter {A : Type}
|
|
theorem T2 ⦃a b : A⦄ (H : a = b) : b = a
|
|
:= symm H
|
|
parameters x y : A
|
|
hypothesis H : x = y
|
|
check T2 H
|
|
check T2
|
|
end
|