src/HOL/ex/Coercion_Examples.thy
changeset 67399 eab6ce8368fa
parent 55932 68c5104d2204
--- a/src/HOL/ex/Coercion_Examples.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/ex/Coercion_Examples.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -65,7 +65,7 @@
 
 term "(1::nat) = (True = (1::nat))"
 
-term "op = (True = (1::nat))"
+term "(=) (True = (1::nat))"
 
 term "[1::nat,True]"