src/HOL/ex/mesontest2.thy
author paulson
Sat, 10 Feb 2007 16:43:23 +0100
changeset 22307 bb31094b4879
parent 19668 6afaf300cb78
child 23774 07968f8cc662
permissions -rw-r--r--
Completing the bug fix from the previous update: the result of unifying type variables must be normalized WRT itself; otherwise instantiation is wrong

(*ID:         $Id$*)
header {* Meson test cases *}

theory mesontest2 imports Main begin

hide const subset

end