src/HOL/Nitpick_Examples/Core_Nits.thy
changeset 67613 ce654b0e6d69
parent 67399 eab6ce8368fa
child 74641 6f801e1073fa
--- a/src/HOL/Nitpick_Examples/Core_Nits.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/Nitpick_Examples/Core_Nits.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -55,7 +55,7 @@
 nitpick [card = 1, expect = genuine]
 oops
 
-lemma "{(a::'a\<times>'a, b::'b)}^-1 = {(b, a)}"
+lemma "{(a::'a\<times>'a, b::'b)}\<inverse> = {(b, a)}"
 nitpick [card = 1-12, expect = none]
 by auto