# HG changeset patch # User wenzelm # Date 1332927974 -7200 # Node ID 6b906beec36ff41143dc2e1ed0eb933d20446ab6 # Parent b9b2e183e94d058a94db24633adbf6577a33ea33 tuned whitespace; diff -r b9b2e183e94d -r 6b906beec36f src/HOL/Unix/Unix.thy --- a/src/HOL/Unix/Unix.thy Wed Mar 28 11:17:32 2012 +0200 +++ b/src/HOL/Unix/Unix.thy Wed Mar 28 11:46:14 2012 +0200 @@ -558,7 +558,7 @@ *} lemma transitions_invariant: - assumes r: "\r x r'. r \x\ r' \ Q r \ P x \ Q r'" + assumes r: "\r x r'. r \x\ r' \ Q r \ P x \ Q r'" and trans: "root =xs\ root'" shows "Q root \ \x \ set xs. P x \ Q root'" using trans